rune/runtime/
function.rs

1use core::fmt;
2use core::future::Future;
3
4use ::rust_alloc::sync::Arc;
5
6use crate as rune;
7use crate::alloc::fmt::TryWrite;
8use crate::alloc::prelude::*;
9use crate::alloc::{self, Box, Vec};
10use crate::function;
11use crate::runtime;
12use crate::runtime::vm::Isolated;
13use crate::shared::AssertSend;
14use crate::Any;
15use crate::Hash;
16
17use super::{
18    Args, Call, ConstValue, Dynamic, Formatter, FromValue, FunctionHandler, GuardedArgs,
19    InstAddress, Output, OwnedTuple, Rtti, RuntimeContext, RuntimeError, Stack, Unit, Value, Vm,
20    VmCall, VmErrorKind, VmHalt, VmResult,
21};
22
23/// The type of a function in Rune.
24///
25/// Functions can be called using call expression syntax, such as `<expr>()`.
26///
27/// There are multiple different kind of things which can be coerced into a
28/// function in Rune:
29/// * Regular functions.
30/// * Closures (which might or might not capture their environment).
31/// * Built-in constructors for tuple types (tuple structs, tuple variants).
32///
33/// # Examples
34///
35/// ```rune
36/// // Captures the constructor for the `Some(<value>)` tuple variant.
37/// let build_some = Some;
38/// assert_eq!(build_some(42), Some(42));
39///
40/// fn build(value) {
41///     Some(value)
42/// }
43///
44/// // Captures the function previously defined.
45/// let build_some = build;
46/// assert_eq!(build_some(42), Some(42));
47/// ```
48#[derive(Any, TryClone)]
49#[repr(transparent)]
50#[rune(item = ::std::ops)]
51pub struct Function(FunctionImpl<Value>);
52
53impl Function {
54    /// Construct a [Function] from a Rust closure.
55    ///
56    /// # Examples
57    ///
58    /// ```
59    /// use rune::{Hash, Vm};
60    /// use rune::runtime::Function;
61    /// use std::sync::Arc;
62    ///
63    /// let mut sources = rune::sources! {
64    ///     entry => {
65    ///         pub fn main(function) {
66    ///             function(41)
67    ///         }
68    ///     }
69    /// };
70    ///
71    /// let unit = rune::prepare(&mut sources).build()?;
72    /// let mut vm = Vm::without_runtime(Arc::new(unit));
73    ///
74    /// let function = Function::new(|value: u32| value + 1);
75    ///
76    /// assert_eq!(function.type_hash(), Hash::EMPTY);
77    ///
78    /// let value = vm.call(["main"], (function,))?;
79    /// let value: u32 = rune::from_value(value)?;
80    /// assert_eq!(value, 42);
81    /// # Ok::<_, rune::support::Error>(())
82    /// ```
83    ///
84    /// Asynchronous functions:
85    ///
86    /// ```
87    /// use rune::{Hash, Vm};
88    /// use rune::runtime::Function;
89    /// use std::sync::Arc;
90    ///
91    /// # futures_executor::block_on(async move {
92    /// let mut sources = rune::sources! {
93    ///     entry => {
94    ///         pub async fn main(function) {
95    ///             function(41).await
96    ///         }
97    ///     }
98    /// };
99    ///
100    /// let unit = rune::prepare(&mut sources).build()?;
101    /// let mut vm = Vm::without_runtime(Arc::new(unit));
102    ///
103    /// let function = Function::new(|value: u32| async move { value + 1 });
104    ///
105    /// assert_eq!(function.type_hash(), Hash::EMPTY);
106    ///
107    /// let value = vm.async_call(["main"], (function,)).await?;
108    /// let value: u32 = rune::from_value(value)?;
109    /// assert_eq!(value, 42);
110    /// # Ok::<_, rune::support::Error>(())
111    /// # })?;
112    /// # Ok::<_, rune::support::Error>(())
113    /// ```
114    pub fn new<F, A, K>(f: F) -> Self
115    where
116        F: function::Function<A, K>,
117        K: function::FunctionKind,
118    {
119        Self(FunctionImpl {
120            inner: Inner::FnHandler(FnHandler {
121                handler: Arc::new(move |stack, addr, args, output| {
122                    f.fn_call(stack, addr, args, output)
123                }),
124                hash: Hash::EMPTY,
125            }),
126        })
127    }
128
129    /// See [`Function::new`].
130    #[deprecated = "Use Function::new() instead"]
131    pub fn function<F, A, K>(f: F) -> Self
132    where
133        F: function::Function<A, K>,
134        K: function::FunctionKind,
135    {
136        Self::new(f)
137    }
138
139    /// See [`Function::function`].
140    #[deprecated = "Use Function::new() instead"]
141    pub fn async_function<F, A>(f: F) -> Self
142    where
143        F: function::Function<A, function::Async>,
144    {
145        Self::new(f)
146    }
147
148    /// Perform an asynchronous call over the function which also implements
149    /// [Send].
150    pub async fn async_send_call<A, T>(&self, args: A) -> VmResult<T>
151    where
152        A: Send + GuardedArgs,
153        T: Send + FromValue,
154    {
155        self.0.async_send_call(args).await
156    }
157
158    /// Perform a call over the function represented by this function pointer.
159    ///
160    /// # Examples
161    ///
162    /// ```
163    /// use rune::{Hash, Vm};
164    /// use rune::runtime::Function;
165    /// use std::sync::Arc;
166    ///
167    /// let mut sources = rune::sources! {
168    ///     entry => {
169    ///         fn add(a, b) {
170    ///             a + b
171    ///         }
172    ///
173    ///         pub fn main() { add }
174    ///     }
175    /// };
176    ///
177    /// let unit = rune::prepare(&mut sources).build()?;
178    /// let mut vm = Vm::without_runtime(Arc::new(unit));
179    /// let value = vm.call(["main"], ())?;
180    ///
181    /// let value: Function = rune::from_value(value)?;
182    /// assert_eq!(value.call::<u32>((1, 2)).into_result()?, 3);
183    /// # Ok::<_, rune::support::Error>(())
184    /// ```
185    pub fn call<T>(&self, args: impl GuardedArgs) -> VmResult<T>
186    where
187        T: FromValue,
188    {
189        self.0.call(args)
190    }
191
192    /// Call with the given virtual machine. This allows for certain
193    /// optimizations, like avoiding the allocation of a new vm state in case
194    /// the call is internal.
195    ///
196    /// A stop reason will be returned in case the function call results in
197    /// a need to suspend the execution.
198    pub(crate) fn call_with_vm(
199        &self,
200        vm: &mut Vm,
201        addr: InstAddress,
202        args: usize,
203        out: Output,
204    ) -> VmResult<Option<VmHalt>> {
205        self.0.call_with_vm(vm, addr, args, out)
206    }
207
208    /// Create a function pointer from a handler.
209    pub(crate) fn from_handler(handler: Arc<FunctionHandler>, hash: Hash) -> Self {
210        Self(FunctionImpl::from_handler(handler, hash))
211    }
212
213    /// Create a function pointer from an offset.
214    pub(crate) fn from_vm_offset(
215        context: Arc<RuntimeContext>,
216        unit: Arc<Unit>,
217        offset: usize,
218        call: Call,
219        args: usize,
220        hash: Hash,
221    ) -> Self {
222        Self(FunctionImpl::from_offset(
223            context, unit, offset, call, args, hash,
224        ))
225    }
226
227    /// Create a function pointer from an offset.
228    pub(crate) fn from_vm_closure(
229        context: Arc<RuntimeContext>,
230        unit: Arc<Unit>,
231        offset: usize,
232        call: Call,
233        args: usize,
234        environment: Box<[Value]>,
235        hash: Hash,
236    ) -> Self {
237        Self(FunctionImpl::from_closure(
238            context,
239            unit,
240            offset,
241            call,
242            args,
243            environment,
244            hash,
245        ))
246    }
247
248    /// Create a function pointer from an offset.
249    pub(crate) fn from_unit_struct(rtti: Arc<Rtti>) -> Self {
250        Self(FunctionImpl::from_unit_struct(rtti))
251    }
252
253    /// Create a function pointer from an offset.
254    pub(crate) fn from_tuple_struct(rtti: Arc<Rtti>, args: usize) -> Self {
255        Self(FunctionImpl::from_tuple_struct(rtti, args))
256    }
257
258    /// Type [Hash][struct@Hash] of the underlying function.
259    ///
260    /// # Examples
261    ///
262    /// The type hash of a top-level function matches what you get out of
263    /// [Hash::type_hash].
264    ///
265    /// ```
266    /// use rune::{Hash, Vm};
267    /// use rune::runtime::Function;
268    /// use std::sync::Arc;
269    ///
270    /// let mut sources = rune::sources! {
271    ///     entry => {
272    ///         fn pony() { }
273    ///
274    ///         pub fn main() { pony }
275    ///     }
276    /// };
277    ///
278    /// let unit = rune::prepare(&mut sources).build()?;
279    /// let mut vm = Vm::without_runtime(Arc::new(unit));
280    /// let pony = vm.call(["main"], ())?;
281    /// let pony: Function = rune::from_value(pony)?;
282    ///
283    /// assert_eq!(pony.type_hash(), Hash::type_hash(["pony"]));
284    /// # Ok::<_, rune::support::Error>(())
285    /// ```
286    pub fn type_hash(&self) -> Hash {
287        self.0.type_hash()
288    }
289
290    /// Try to convert into a [SyncFunction]. This might not be possible if this
291    /// function is something which is not [Sync], like a closure capturing
292    /// context which is not thread-safe.
293    ///
294    /// # Examples
295    ///
296    /// ```
297    /// use rune::{Hash, Vm};
298    /// use rune::runtime::Function;
299    /// use std::sync::Arc;
300    ///
301    /// let mut sources = rune::sources! {
302    ///     entry => {
303    ///         fn pony() { }
304    ///
305    ///         pub fn main() { pony }
306    ///     }
307    /// };
308    ///
309    /// let unit = rune::prepare(&mut sources).build()?;
310    /// let mut vm = Vm::without_runtime(Arc::new(unit));
311    /// let pony = vm.call(["main"], ())?;
312    /// let pony: Function = rune::from_value(pony)?;
313    ///
314    /// // This is fine, since `pony` is a free function.
315    /// let pony = pony.into_sync()?;
316    ///
317    /// assert_eq!(pony.type_hash(), Hash::type_hash(["pony"]));
318    /// # Ok::<_, rune::support::Error>(())
319    /// ```
320    ///
321    /// The following *does not* work, because we return a closure which tries
322    /// to make use of a [Generator][crate::runtime::Generator] which is not a
323    /// constant value.
324    ///
325    /// ```
326    /// use rune::{Hash, Vm};
327    /// use rune::runtime::Function;
328    /// use std::sync::Arc;
329    ///
330    /// let mut sources = rune::sources! {
331    ///     entry => {
332    ///         fn generator() {
333    ///             yield 42;
334    ///         }
335    ///
336    ///         pub fn main() {
337    ///             let g = generator();
338    ///
339    ///             move || {
340    ///                 g.next()
341    ///             }
342    ///         }
343    ///     }
344    /// };
345    ///
346    /// let unit = rune::prepare(&mut sources).build()?;
347    /// let mut vm = Vm::without_runtime(Arc::new(unit));
348    /// let closure = vm.call(["main"], ())?;
349    /// let closure: Function = rune::from_value(closure)?;
350    ///
351    /// // This is *not* fine since the returned closure has captured a
352    /// // generator which is not a constant value.
353    /// assert!(closure.into_sync().is_err());
354    /// # Ok::<_, rune::support::Error>(())
355    /// ```
356    pub fn into_sync(self) -> Result<SyncFunction, RuntimeError> {
357        Ok(SyncFunction(self.0.into_sync()?))
358    }
359
360    /// Clone a function.
361    ///
362    /// # Examples
363    ///
364    /// ```rune
365    /// fn function() {
366    ///     42
367    /// }
368    ///
369    /// let a = function;
370    /// let b = a.clone();
371    /// assert_eq!(a(), b());
372    /// ```
373    #[rune::function(keep, protocol = CLONE)]
374    fn clone(&self) -> VmResult<Function> {
375        VmResult::Ok(vm_try!(self.try_clone()))
376    }
377
378    /// Debug format a function.
379    ///
380    /// # Examples
381    ///
382    /// ```rune
383    /// fn function() {
384    ///     42
385    /// }
386    ///
387    /// println!("{function:?}");
388    /// ``
389    #[rune::function(keep, protocol = DEBUG_FMT)]
390    fn debug_fmt(&self, f: &mut Formatter) -> VmResult<()> {
391        vm_write!(f, "{self:?}")
392    }
393}
394
395/// A callable sync function. This currently only supports a subset of values
396/// that are supported by the Vm.
397#[repr(transparent)]
398pub struct SyncFunction(FunctionImpl<ConstValue>);
399
400assert_impl!(SyncFunction: Send + Sync);
401
402impl SyncFunction {
403    /// Perform an asynchronous call over the function which also implements
404    /// [Send].
405    ///
406    /// # Examples
407    ///
408    /// ```
409    /// use rune::{Hash, Vm};
410    /// use rune::runtime::SyncFunction;
411    /// use std::sync::Arc;
412    ///
413    /// # futures_executor::block_on(async move {
414    /// let mut sources = rune::sources! {
415    ///     entry => {
416    ///         async fn add(a, b) {
417    ///             a + b
418    ///         }
419    ///
420    ///         pub fn main() { add }
421    ///     }
422    /// };
423    ///
424    /// let unit = rune::prepare(&mut sources).build()?;
425    /// let mut vm = Vm::without_runtime(Arc::new(unit));
426    /// let add = vm.call(["main"], ())?;
427    /// let add: SyncFunction = rune::from_value(add)?;
428    ///
429    /// let value = add.async_send_call::<u32>((1, 2)).await.into_result()?;
430    /// assert_eq!(value, 3);
431    /// # Ok::<_, rune::support::Error>(())
432    /// # })?;
433    /// # Ok::<_, rune::support::Error>(())
434    /// ```
435    pub async fn async_send_call<T>(&self, args: impl GuardedArgs + Send) -> VmResult<T>
436    where
437        T: Send + FromValue,
438    {
439        self.0.async_send_call(args).await
440    }
441
442    /// Perform a call over the function represented by this function pointer.
443    ///
444    /// # Examples
445    ///
446    /// ```
447    /// use rune::{Hash, Vm};
448    /// use rune::runtime::SyncFunction;
449    /// use std::sync::Arc;
450    ///
451    /// let mut sources = rune::sources! {
452    ///     entry => {
453    ///         fn add(a, b) {
454    ///             a + b
455    ///         }
456    ///
457    ///         pub fn main() { add }
458    ///     }
459    /// };
460    ///
461    /// let unit = rune::prepare(&mut sources).build()?;
462    /// let mut vm = Vm::without_runtime(Arc::new(unit));
463    /// let add = vm.call(["main"], ())?;
464    /// let add: SyncFunction = rune::from_value(add)?;
465    ///
466    /// assert_eq!(add.call::<u32>((1, 2)).into_result()?, 3);
467    /// # Ok::<_, rune::support::Error>(())
468    /// ```
469    pub fn call<T>(&self, args: impl GuardedArgs) -> VmResult<T>
470    where
471        T: FromValue,
472    {
473        self.0.call(args)
474    }
475
476    /// Type [Hash][struct@Hash] of the underlying function.
477    ///
478    /// # Examples
479    ///
480    /// The type hash of a top-level function matches what you get out of
481    /// [Hash::type_hash].
482    ///
483    /// ```
484    /// use rune::{Hash, Vm};
485    /// use rune::runtime::SyncFunction;
486    /// use std::sync::Arc;
487    ///
488    /// let mut sources = rune::sources! {
489    ///     entry => {
490    ///         fn pony() { }
491    ///
492    ///         pub fn main() { pony }
493    ///     }
494    /// };
495    ///
496    /// let unit = rune::prepare(&mut sources).build()?;
497    /// let mut vm = Vm::without_runtime(Arc::new(unit));
498    /// let pony = vm.call(["main"], ())?;
499    /// let pony: SyncFunction = rune::from_value(pony)?;
500    ///
501    /// assert_eq!(pony.type_hash(), Hash::type_hash(["pony"]));
502    /// # Ok::<_, rune::support::Error>(())
503    /// ```
504    pub fn type_hash(&self) -> Hash {
505        self.0.type_hash()
506    }
507}
508
509impl TryClone for SyncFunction {
510    fn try_clone(&self) -> alloc::Result<Self> {
511        Ok(Self(self.0.try_clone()?))
512    }
513}
514
515/// A stored function, of some specific kind.
516struct FunctionImpl<V> {
517    inner: Inner<V>,
518}
519
520impl<V> TryClone for FunctionImpl<V>
521where
522    V: TryClone,
523{
524    #[inline]
525    fn try_clone(&self) -> alloc::Result<Self> {
526        Ok(Self {
527            inner: self.inner.try_clone()?,
528        })
529    }
530}
531
532impl<V> FunctionImpl<V>
533where
534    V: TryClone,
535    OwnedTuple: TryFrom<Box<[V]>>,
536    VmErrorKind: From<<OwnedTuple as TryFrom<Box<[V]>>>::Error>,
537{
538    fn call<T>(&self, args: impl GuardedArgs) -> VmResult<T>
539    where
540        T: FromValue,
541    {
542        let value = match &self.inner {
543            Inner::FnHandler(handler) => {
544                let count = args.count();
545                let size = count.max(1);
546                // Ensure we have space for the return value.
547                let mut stack = vm_try!(Stack::with_capacity(size));
548                let _guard = vm_try!(unsafe { args.guarded_into_stack(&mut stack) });
549                vm_try!(stack.resize(size));
550                vm_try!((handler.handler)(
551                    &mut stack,
552                    InstAddress::ZERO,
553                    count,
554                    InstAddress::ZERO.output()
555                ));
556                stack.at(InstAddress::ZERO).clone()
557            }
558            Inner::FnOffset(fn_offset) => {
559                vm_try!(fn_offset.call(args, ()))
560            }
561            Inner::FnClosureOffset(closure) => {
562                let environment = vm_try!(closure.environment.try_clone());
563                let environment = vm_try!(OwnedTuple::try_from(environment));
564                vm_try!(closure.fn_offset.call(args, (environment,)))
565            }
566            Inner::FnUnitStruct(empty) => {
567                vm_try!(check_args(args.count(), 0));
568                vm_try!(Value::empty_struct(empty.rtti.clone()))
569            }
570            Inner::FnTupleStruct(tuple) => {
571                vm_try!(check_args(args.count(), tuple.args));
572                // SAFETY: We don't let the guard outlive the value.
573                let (args, _guard) = vm_try!(unsafe { args.guarded_into_vec() });
574                vm_try!(Value::tuple_struct(tuple.rtti.clone(), args))
575            }
576        };
577
578        VmResult::Ok(vm_try!(T::from_value(value)))
579    }
580
581    fn async_send_call<'a, A, T>(&'a self, args: A) -> impl Future<Output = VmResult<T>> + Send + 'a
582    where
583        A: 'a + Send + GuardedArgs,
584        T: 'a + Send + FromValue,
585    {
586        let future = async move {
587            let value: Value = vm_try!(self.call(args));
588
589            let value = match vm_try!(value.try_borrow_mut::<runtime::Future>()) {
590                Some(future) => vm_try!(future.await),
591                None => value,
592            };
593
594            VmResult::Ok(vm_try!(T::from_value(value)))
595        };
596
597        // Safety: Future is send because there is no way to call this
598        // function in a manner which allows any values from the future
599        // to escape outside of this future, hence it can only be
600        // scheduled by one thread at a time.
601        unsafe { AssertSend::new(future) }
602    }
603
604    /// Call with the given virtual machine. This allows for certain
605    /// optimizations, like avoiding the allocation of a new vm state in case
606    /// the call is internal.
607    ///
608    /// A stop reason will be returned in case the function call results in
609    /// a need to suspend the execution.
610    pub(crate) fn call_with_vm(
611        &self,
612        vm: &mut Vm,
613        addr: InstAddress,
614        args: usize,
615        out: Output,
616    ) -> VmResult<Option<VmHalt>> {
617        let reason = match &self.inner {
618            Inner::FnHandler(handler) => {
619                vm_try!((handler.handler)(vm.stack_mut(), addr, args, out));
620                None
621            }
622            Inner::FnOffset(fn_offset) => {
623                if let Some(vm_call) = vm_try!(fn_offset.call_with_vm(vm, addr, args, (), out)) {
624                    return VmResult::Ok(Some(VmHalt::VmCall(vm_call)));
625                }
626
627                None
628            }
629            Inner::FnClosureOffset(closure) => {
630                let environment = vm_try!(closure.environment.try_clone());
631                let environment = vm_try!(OwnedTuple::try_from(environment));
632
633                if let Some(vm_call) =
634                    vm_try!(closure
635                        .fn_offset
636                        .call_with_vm(vm, addr, args, (environment,), out))
637                {
638                    return VmResult::Ok(Some(VmHalt::VmCall(vm_call)));
639                }
640
641                None
642            }
643            Inner::FnUnitStruct(empty) => {
644                vm_try!(check_args(args, 0));
645                vm_try!(out.store(vm.stack_mut(), || Value::empty_struct(empty.rtti.clone())));
646                None
647            }
648            Inner::FnTupleStruct(tuple) => {
649                vm_try!(check_args(args, tuple.args));
650
651                let seq = vm_try!(vm.stack().slice_at(addr, args));
652                let data = seq.iter().cloned();
653                let value = vm_try!(Dynamic::new(tuple.rtti.clone(), data));
654                vm_try!(out.store(vm.stack_mut(), value));
655                None
656            }
657        };
658
659        VmResult::Ok(reason)
660    }
661
662    /// Create a function pointer from a handler.
663    pub(crate) fn from_handler(handler: Arc<FunctionHandler>, hash: Hash) -> Self {
664        Self {
665            inner: Inner::FnHandler(FnHandler { handler, hash }),
666        }
667    }
668
669    /// Create a function pointer from an offset.
670    pub(crate) fn from_offset(
671        context: Arc<RuntimeContext>,
672        unit: Arc<Unit>,
673        offset: usize,
674        call: Call,
675        args: usize,
676        hash: Hash,
677    ) -> Self {
678        Self {
679            inner: Inner::FnOffset(FnOffset {
680                context,
681                unit,
682                offset,
683                call,
684                args,
685                hash,
686            }),
687        }
688    }
689
690    /// Create a function pointer from an offset.
691    pub(crate) fn from_closure(
692        context: Arc<RuntimeContext>,
693        unit: Arc<Unit>,
694        offset: usize,
695        call: Call,
696        args: usize,
697        environment: Box<[V]>,
698        hash: Hash,
699    ) -> Self {
700        Self {
701            inner: Inner::FnClosureOffset(FnClosureOffset {
702                fn_offset: FnOffset {
703                    context,
704                    unit,
705                    offset,
706                    call,
707                    args,
708                    hash,
709                },
710                environment,
711            }),
712        }
713    }
714
715    /// Create a function pointer from an offset.
716    pub(crate) fn from_unit_struct(rtti: Arc<Rtti>) -> Self {
717        Self {
718            inner: Inner::FnUnitStruct(FnUnitStruct { rtti }),
719        }
720    }
721
722    /// Create a function pointer from an offset.
723    pub(crate) fn from_tuple_struct(rtti: Arc<Rtti>, args: usize) -> Self {
724        Self {
725            inner: Inner::FnTupleStruct(FnTupleStruct { rtti, args }),
726        }
727    }
728
729    #[inline]
730    fn type_hash(&self) -> Hash {
731        match &self.inner {
732            Inner::FnHandler(FnHandler { hash, .. }) | Inner::FnOffset(FnOffset { hash, .. }) => {
733                *hash
734            }
735            Inner::FnClosureOffset(fco) => fco.fn_offset.hash,
736            Inner::FnUnitStruct(func) => func.rtti.type_hash(),
737            Inner::FnTupleStruct(func) => func.rtti.type_hash(),
738        }
739    }
740}
741
742impl FunctionImpl<Value> {
743    /// Try to convert into a [SyncFunction].
744    fn into_sync(self) -> Result<FunctionImpl<ConstValue>, RuntimeError> {
745        let inner = match self.inner {
746            Inner::FnClosureOffset(closure) => {
747                let mut env = Vec::try_with_capacity(closure.environment.len())?;
748
749                for value in Vec::from(closure.environment) {
750                    env.try_push(FromValue::from_value(value)?)?;
751                }
752
753                Inner::FnClosureOffset(FnClosureOffset {
754                    fn_offset: closure.fn_offset,
755                    environment: env.try_into_boxed_slice()?,
756                })
757            }
758            Inner::FnHandler(inner) => Inner::FnHandler(inner),
759            Inner::FnOffset(inner) => Inner::FnOffset(inner),
760            Inner::FnUnitStruct(inner) => Inner::FnUnitStruct(inner),
761            Inner::FnTupleStruct(inner) => Inner::FnTupleStruct(inner),
762        };
763
764        Ok(FunctionImpl { inner })
765    }
766}
767
768impl fmt::Debug for Function {
769    fn fmt(&self, f: &mut fmt::Formatter<'_>) -> fmt::Result {
770        match &self.0.inner {
771            Inner::FnHandler(handler) => {
772                write!(f, "native function ({:p})", handler.handler.as_ref())?;
773            }
774            Inner::FnOffset(offset) => {
775                write!(f, "{} function (at: 0x{:x})", offset.call, offset.offset)?;
776            }
777            Inner::FnClosureOffset(closure) => {
778                write!(
779                    f,
780                    "closure (at: 0x{:x}, env:{:?})",
781                    closure.fn_offset.offset, closure.environment
782                )?;
783            }
784            Inner::FnUnitStruct(empty) => {
785                write!(f, "empty {}", empty.rtti.item)?;
786            }
787            Inner::FnTupleStruct(tuple) => {
788                write!(f, "tuple {}", tuple.rtti.item)?;
789            }
790        }
791
792        Ok(())
793    }
794}
795
796#[derive(Debug)]
797enum Inner<V> {
798    /// A native function handler.
799    /// This is wrapped as an `Arc<dyn FunctionHandler>`.
800    FnHandler(FnHandler),
801    /// The offset to a free function.
802    ///
803    /// This also captures the context and unit it belongs to allow for external
804    /// calls.
805    FnOffset(FnOffset),
806    /// A closure with a captured environment.
807    ///
808    /// This also captures the context and unit it belongs to allow for external
809    /// calls.
810    FnClosureOffset(FnClosureOffset<V>),
811    /// Constructor for a unit struct.
812    FnUnitStruct(FnUnitStruct),
813    /// Constructor for a tuple.
814    FnTupleStruct(FnTupleStruct),
815}
816
817impl<V> TryClone for Inner<V>
818where
819    V: TryClone,
820{
821    fn try_clone(&self) -> alloc::Result<Self> {
822        Ok(match self {
823            Inner::FnHandler(inner) => Inner::FnHandler(inner.clone()),
824            Inner::FnOffset(inner) => Inner::FnOffset(inner.clone()),
825            Inner::FnClosureOffset(inner) => Inner::FnClosureOffset(inner.try_clone()?),
826            Inner::FnUnitStruct(inner) => Inner::FnUnitStruct(inner.clone()),
827            Inner::FnTupleStruct(inner) => Inner::FnTupleStruct(inner.clone()),
828        })
829    }
830}
831
832#[derive(Clone, TryClone)]
833struct FnHandler {
834    /// The function handler.
835    handler: Arc<FunctionHandler>,
836    /// Hash for the function type
837    hash: Hash,
838}
839
840impl fmt::Debug for FnHandler {
841    fn fmt(&self, f: &mut fmt::Formatter<'_>) -> fmt::Result {
842        write!(f, "FnHandler")
843    }
844}
845
846#[derive(Clone, TryClone)]
847struct FnOffset {
848    context: Arc<RuntimeContext>,
849    /// The unit where the function resides.
850    unit: Arc<Unit>,
851    /// The offset of the function.
852    offset: usize,
853    /// The calling convention.
854    call: Call,
855    /// The number of arguments the function takes.
856    args: usize,
857    /// Hash for the function type
858    hash: Hash,
859}
860
861impl FnOffset {
862    /// Perform a call into the specified offset and return the produced value.
863    #[tracing::instrument(skip_all, fields(args = args.count(), extra = extra.count(), ?self.offset, ?self.call, ?self.args, ?self.hash))]
864    fn call(&self, args: impl GuardedArgs, extra: impl Args) -> VmResult<Value> {
865        vm_try!(check_args(
866            args.count().wrapping_add(extra.count()),
867            self.args
868        ));
869
870        let mut vm = Vm::new(self.context.clone(), self.unit.clone());
871
872        vm.set_ip(self.offset);
873        let _guard = vm_try!(unsafe { args.guarded_into_stack(vm.stack_mut()) });
874        vm_try!(extra.into_stack(vm.stack_mut()));
875
876        self.call.call_with_vm(vm)
877    }
878
879    /// Perform a potentially optimized call into the specified vm.
880    ///
881    /// This will cause a halt in case the vm being called into isn't the same
882    /// as the context and unit of the function.
883    #[tracing::instrument(skip_all, fields(args, extra = extra.count(), keep, ?self.offset, ?self.call, ?self.args, ?self.hash))]
884    fn call_with_vm(
885        &self,
886        vm: &mut Vm,
887        addr: InstAddress,
888        args: usize,
889        extra: impl Args,
890        out: Output,
891    ) -> VmResult<Option<VmCall>> {
892        vm_try!(check_args(args.wrapping_add(extra.count()), self.args));
893
894        let same_unit = matches!(self.call, Call::Immediate if vm.is_same_unit(&self.unit));
895        let same_context =
896            matches!(self.call, Call::Immediate if vm.is_same_context(&self.context));
897
898        vm_try!(vm.push_call_frame(self.offset, addr, args, Isolated::new(!same_context), out));
899        vm_try!(extra.into_stack(vm.stack_mut()));
900
901        // Fast path, just allocate a call frame and keep running.
902        if same_context && same_unit {
903            tracing::trace!("same context and unit");
904            return VmResult::Ok(None);
905        }
906
907        VmResult::Ok(Some(VmCall::new(
908            self.call,
909            (!same_context).then(|| self.context.clone()),
910            (!same_unit).then(|| self.unit.clone()),
911            out,
912        )))
913    }
914}
915
916impl fmt::Debug for FnOffset {
917    fn fmt(&self, f: &mut fmt::Formatter<'_>) -> fmt::Result {
918        f.debug_struct("FnOffset")
919            .field("context", &(&self.context as *const _))
920            .field("unit", &(&self.unit as *const _))
921            .field("offset", &self.offset)
922            .field("call", &self.call)
923            .field("args", &self.args)
924            .finish()
925    }
926}
927
928#[derive(Debug)]
929struct FnClosureOffset<V> {
930    /// The offset in the associated unit that the function lives.
931    fn_offset: FnOffset,
932    /// Captured environment.
933    environment: Box<[V]>,
934}
935
936impl<V> TryClone for FnClosureOffset<V>
937where
938    V: TryClone,
939{
940    #[inline]
941    fn try_clone(&self) -> alloc::Result<Self> {
942        Ok(Self {
943            fn_offset: self.fn_offset.clone(),
944            environment: self.environment.try_clone()?,
945        })
946    }
947}
948
949#[derive(Debug, Clone, TryClone)]
950struct FnUnitStruct {
951    /// The type of the empty.
952    rtti: Arc<Rtti>,
953}
954
955#[derive(Debug, Clone, TryClone)]
956struct FnTupleStruct {
957    /// The type of the tuple.
958    rtti: Arc<Rtti>,
959    /// The number of arguments the tuple takes.
960    args: usize,
961}
962
963impl FromValue for SyncFunction {
964    #[inline]
965    fn from_value(value: Value) -> Result<Self, RuntimeError> {
966        value.downcast::<Function>()?.into_sync()
967    }
968}
969
970fn check_args(actual: usize, expected: usize) -> VmResult<()> {
971    if actual != expected {
972        return VmResult::err(VmErrorKind::BadArgumentCount { expected, actual });
973    }
974
975    VmResult::Ok(())
976}