summaryrefslogtreecommitdiff
path: root/tests/lean/Traits.lean
diff options
context:
space:
mode:
authorSon Ho2023-11-21 14:57:38 +0100
committerSon Ho2023-11-21 14:57:38 +0100
commit137cc7335e64fcb70c254e7fd2a6fa353fb43e61 (patch)
treef703dc52640670ad9e634ea0d6cc93c0c98cbede /tests/lean/Traits.lean
parentd564a010893653edea0df518e0b740fadf7df031 (diff)
Regenerate the files
Diffstat (limited to 'tests/lean/Traits.lean')
-rw-r--r--tests/lean/Traits.lean219
1 files changed, 146 insertions, 73 deletions
diff --git a/tests/lean/Traits.lean b/tests/lean/Traits.lean
index 51a05581..f854da76 100644
--- a/tests/lean/Traits.lean
+++ b/tests/lean/Traits.lean
@@ -5,25 +5,30 @@ open Primitives
namespace traits
-/- Trait declaration: [traits::BoolTrait] -/
+/- Trait declaration: [traits::BoolTrait]
+ Source: 'src/traits.rs', lines 1:0-1:19 -/
structure BoolTrait (Self : Type) where
get_bool : Self → Result Bool
-/- [traits::{bool}::get_bool]: forward function -/
+/- [traits::{bool}::get_bool]: forward function
+ Source: 'src/traits.rs', lines 12:4-12:30 -/
def Bool.get_bool (self : Bool) : Result Bool :=
Result.ret self
-/- Trait implementation: [traits::{bool}] -/
+/- Trait implementation: [traits::{bool}]
+ Source: 'src/traits.rs', lines 11:0-11:23 -/
def traits.BoolTraitBoolInst : BoolTrait Bool := {
get_bool := Bool.get_bool
}
-/- [traits::BoolTrait::ret_true]: forward function -/
+/- [traits::BoolTrait::ret_true]: forward function
+ Source: 'src/traits.rs', lines 6:4-6:30 -/
def BoolTrait.ret_true
{Self : Type} (self_clause : BoolTrait Self) (self : Self) : Result Bool :=
Result.ret true
-/- [traits::test_bool_trait_bool]: forward function -/
+/- [traits::test_bool_trait_bool]: forward function
+ Source: 'src/traits.rs', lines 17:0-17:44 -/
def test_bool_trait_bool (x : Bool) : Result Bool :=
do
let b ← Bool.get_bool x
@@ -31,19 +36,22 @@ def test_bool_trait_bool (x : Bool) : Result Bool :=
then BoolTrait.ret_true traits.BoolTraitBoolInst x
else Result.ret false
-/- [traits::{core::option::Option<T>#1}::get_bool]: forward function -/
+/- [traits::{core::option::Option<T>#1}::get_bool]: forward function
+ Source: 'src/traits.rs', lines 23:4-23:30 -/
def Option.get_bool (T : Type) (self : Option T) : Result Bool :=
match self with
| none => Result.ret false
| some t => Result.ret true
-/- Trait implementation: [traits::{core::option::Option<T>#1}] -/
+/- Trait implementation: [traits::{core::option::Option<T>#1}]
+ Source: 'src/traits.rs', lines 22:0-22:31 -/
def traits.BoolTraitcoreoptionOptionTInst (T : Type) : BoolTrait (Option T)
:= {
get_bool := Option.get_bool T
}
-/- [traits::test_bool_trait_option]: forward function -/
+/- [traits::test_bool_trait_option]: forward function
+ Source: 'src/traits.rs', lines 31:0-31:54 -/
def test_bool_trait_option (T : Type) (x : Option T) : Result Bool :=
do
let b ← Option.get_bool T x
@@ -51,24 +59,29 @@ def test_bool_trait_option (T : Type) (x : Option T) : Result Bool :=
then BoolTrait.ret_true (traits.BoolTraitcoreoptionOptionTInst T) x
else Result.ret false
-/- [traits::test_bool_trait]: forward function -/
+/- [traits::test_bool_trait]: forward function
+ Source: 'src/traits.rs', lines 35:0-35:50 -/
def test_bool_trait (T : Type) (inst : BoolTrait T) (x : T) : Result Bool :=
inst.get_bool x
-/- Trait declaration: [traits::ToU64] -/
+/- Trait declaration: [traits::ToU64]
+ Source: 'src/traits.rs', lines 39:0-39:15 -/
structure ToU64 (Self : Type) where
to_u64 : Self → Result U64
-/- [traits::{u64#2}::to_u64]: forward function -/
+/- [traits::{u64#2}::to_u64]: forward function
+ Source: 'src/traits.rs', lines 44:4-44:26 -/
def U64.to_u64 (self : U64) : Result U64 :=
Result.ret self
-/- Trait implementation: [traits::{u64#2}] -/
+/- Trait implementation: [traits::{u64#2}]
+ Source: 'src/traits.rs', lines 43:0-43:18 -/
def traits.ToU64U64Inst : ToU64 U64 := {
to_u64 := U64.to_u64
}
-/- [traits::{(A, A)#3}::to_u64]: forward function -/
+/- [traits::{(A, A)#3}::to_u64]: forward function
+ Source: 'src/traits.rs', lines 50:4-50:26 -/
def Pair.to_u64 (A : Type) (inst : ToU64 A) (self : (A × A)) : Result U64 :=
do
let (t, t0) := self
@@ -76,106 +89,128 @@ def Pair.to_u64 (A : Type) (inst : ToU64 A) (self : (A × A)) : Result U64 :=
let i0 ← inst.to_u64 t0
i + i0
-/- Trait implementation: [traits::{(A, A)#3}] -/
+/- Trait implementation: [traits::{(A, A)#3}]
+ Source: 'src/traits.rs', lines 49:0-49:31 -/
def traits.ToU64TupleAAInst (A : Type) (inst : ToU64 A) : ToU64 (A × A) := {
to_u64 := Pair.to_u64 A inst
}
-/- [traits::f]: forward function -/
+/- [traits::f]: forward function
+ Source: 'src/traits.rs', lines 55:0-55:36 -/
def f (T : Type) (inst : ToU64 T) (x : (T × T)) : Result U64 :=
Pair.to_u64 T inst x
-/- [traits::g]: forward function -/
+/- [traits::g]: forward function
+ Source: 'src/traits.rs', lines 59:0-61:18 -/
def g (T : Type) (inst : ToU64 (T × T)) (x : (T × T)) : Result U64 :=
inst.to_u64 x
-/- [traits::h0]: forward function -/
+/- [traits::h0]: forward function
+ Source: 'src/traits.rs', lines 66:0-66:24 -/
def h0 (x : U64) : Result U64 :=
U64.to_u64 x
-/- [traits::Wrapper] -/
+/- [traits::Wrapper]
+ Source: 'src/traits.rs', lines 70:0-70:21 -/
structure Wrapper (T : Type) where
x : T
-/- [traits::{traits::Wrapper<T>#4}::to_u64]: forward function -/
+/- [traits::{traits::Wrapper<T>#4}::to_u64]: forward function
+ Source: 'src/traits.rs', lines 75:4-75:26 -/
def Wrapper.to_u64
(T : Type) (inst : ToU64 T) (self : Wrapper T) : Result U64 :=
inst.to_u64 self.x
-/- Trait implementation: [traits::{traits::Wrapper<T>#4}] -/
+/- Trait implementation: [traits::{traits::Wrapper<T>#4}]
+ Source: 'src/traits.rs', lines 74:0-74:35 -/
def traits.ToU64traitsWrapperTInst (T : Type) (inst : ToU64 T) : ToU64 (Wrapper
T) := {
to_u64 := Wrapper.to_u64 T inst
}
-/- [traits::h1]: forward function -/
+/- [traits::h1]: forward function
+ Source: 'src/traits.rs', lines 80:0-80:33 -/
def h1 (x : Wrapper U64) : Result U64 :=
Wrapper.to_u64 U64 traits.ToU64U64Inst x
-/- [traits::h2]: forward function -/
+/- [traits::h2]: forward function
+ Source: 'src/traits.rs', lines 84:0-84:41 -/
def h2 (T : Type) (inst : ToU64 T) (x : Wrapper T) : Result U64 :=
Wrapper.to_u64 T inst x
-/- Trait declaration: [traits::ToType] -/
+/- Trait declaration: [traits::ToType]
+ Source: 'src/traits.rs', lines 88:0-88:19 -/
structure ToType (Self T : Type) where
to_type : Self → Result T
-/- [traits::{u64#5}::to_type]: forward function -/
+/- [traits::{u64#5}::to_type]: forward function
+ Source: 'src/traits.rs', lines 93:4-93:28 -/
def U64.to_type (self : U64) : Result Bool :=
Result.ret (self > 0#u64)
-/- Trait implementation: [traits::{u64#5}] -/
+/- Trait implementation: [traits::{u64#5}]
+ Source: 'src/traits.rs', lines 92:0-92:25 -/
def traits.ToTypeU64BoolInst : ToType U64 Bool := {
to_type := U64.to_type
}
-/- Trait declaration: [traits::OfType] -/
+/- Trait declaration: [traits::OfType]
+ Source: 'src/traits.rs', lines 98:0-98:16 -/
structure OfType (Self : Type) where
of_type : forall (T : Type) (inst : ToType T Self), T → Result Self
-/- [traits::h3]: forward function -/
+/- [traits::h3]: forward function
+ Source: 'src/traits.rs', lines 104:0-104:50 -/
def h3
(T1 T2 : Type) (inst : OfType T1) (inst0 : ToType T2 T1) (y : T2) :
Result T1
:=
inst.of_type T2 inst0 y
-/- Trait declaration: [traits::OfTypeBis] -/
+/- Trait declaration: [traits::OfTypeBis]
+ Source: 'src/traits.rs', lines 109:0-109:36 -/
structure OfTypeBis (Self T : Type) where
parent_clause_0 : ToType T Self
of_type : T → Result Self
-/- [traits::h4]: forward function -/
+/- [traits::h4]: forward function
+ Source: 'src/traits.rs', lines 118:0-118:57 -/
def h4
(T1 T2 : Type) (inst : OfTypeBis T1 T2) (inst0 : ToType T2 T1) (y : T2) :
Result T1
:=
inst.of_type y
-/- [traits::TestType] -/
+/- [traits::TestType]
+ Source: 'src/traits.rs', lines 122:0-122:22 -/
structure TestType (T : Type) where
_0 : T
-/- [traits::{traits::TestType<T>#6}::test::TestType1] -/
+/- [traits::{traits::TestType<T>#6}::test::TestType1]
+ Source: 'src/traits.rs', lines 127:8-127:24 -/
structure TestType.test.TestType1 where
_0 : U64
-/- Trait declaration: [traits::{traits::TestType<T>#6}::test::TestTrait] -/
+/- Trait declaration: [traits::{traits::TestType<T>#6}::test::TestTrait]
+ Source: 'src/traits.rs', lines 128:8-128:23 -/
structure TestType.test.TestTrait (Self : Type) where
test : Self → Result Bool
-/- [traits::{traits::TestType<T>#6}::test::{traits::{traits::TestType<T>#6}::test::TestType1}::test]: forward function -/
+/- [traits::{traits::TestType<T>#6}::test::{traits::{traits::TestType<T>#6}::test::TestType1}::test]: forward function
+ Source: 'src/traits.rs', lines 139:12-139:34 -/
def TestType.test.TestType1.test
(self : TestType.test.TestType1) : Result Bool :=
Result.ret (self._0 > 1#u64)
-/- Trait implementation: [traits::{traits::TestType<T>#6}::test::{traits::{traits::TestType<T>#6}::test::TestType1}] -/
+/- Trait implementation: [traits::{traits::TestType<T>#6}::test::{traits::{traits::TestType<T>#6}::test::TestType1}]
+ Source: 'src/traits.rs', lines 138:8-138:36 -/
def traits.TestType.test.TestTraittraitstraitsTestTypeTtestTestType1Inst :
TestType.test.TestTrait TestType.test.TestType1 := {
test := TestType.test.TestType1.test
}
-/- [traits::{traits::TestType<T>#6}::test]: forward function -/
+/- [traits::{traits::TestType<T>#6}::test]: forward function
+ Source: 'src/traits.rs', lines 126:4-126:36 -/
def TestType.test
(T : Type) (inst : ToU64 T) (self : TestType T) (x : T) : Result Bool :=
do
@@ -184,27 +219,32 @@ def TestType.test
then TestType.test.TestType1.test { _0 := 0#u64 }
else Result.ret false
-/- [traits::BoolWrapper] -/
+/- [traits::BoolWrapper]
+ Source: 'src/traits.rs', lines 150:0-150:22 -/
structure BoolWrapper where
_0 : Bool
-/- [traits::{traits::BoolWrapper#7}::to_type]: forward function -/
+/- [traits::{traits::BoolWrapper#7}::to_type]: forward function
+ Source: 'src/traits.rs', lines 156:4-156:25 -/
def BoolWrapper.to_type
(T : Type) (inst : ToType Bool T) (self : BoolWrapper) : Result T :=
inst.to_type self._0
-/- Trait implementation: [traits::{traits::BoolWrapper#7}] -/
+/- Trait implementation: [traits::{traits::BoolWrapper#7}]
+ Source: 'src/traits.rs', lines 152:0-152:33 -/
def traits.ToTypetraitsBoolWrapperTInst (T : Type) (inst : ToType Bool T) :
ToType BoolWrapper T := {
to_type := BoolWrapper.to_type T inst
}
-/- [traits::WithConstTy::LEN2] -/
+/- [traits::WithConstTy::LEN2]
+ Source: 'src/traits.rs', lines 164:4-164:21 -/
def with_const_ty_len2_body : Result Usize := Result.ret 32#usize
def with_const_ty_len2_c : Usize :=
eval_global with_const_ty_len2_body (by simp)
-/- Trait declaration: [traits::WithConstTy] -/
+/- Trait declaration: [traits::WithConstTy]
+ Source: 'src/traits.rs', lines 161:0-161:39 -/
structure WithConstTy (Self : Type) (LEN : Usize) where
LEN1 : Usize
LEN2 : Usize
@@ -213,16 +253,19 @@ structure WithConstTy (Self : Type) (LEN : Usize) where
W_clause_0 : ToU64 W
f : W → Array U8 LEN → Result W
-/- [traits::{bool#8}::LEN1] -/
+/- [traits::{bool#8}::LEN1]
+ Source: 'src/traits.rs', lines 175:4-175:21 -/
def bool_len1_body : Result Usize := Result.ret 12#usize
def bool_len1_c : Usize := eval_global bool_len1_body (by simp)
/- [traits::{bool#8}::f]: merged forward/backward function
- (there is a single backward function, and the forward function returns ()) -/
+ (there is a single backward function, and the forward function returns ())
+ Source: 'src/traits.rs', lines 180:4-180:39 -/
def Bool.f (i : U64) (a : Array U8 32#usize) : Result U64 :=
Result.ret i
-/- Trait implementation: [traits::{bool#8}] -/
+/- Trait implementation: [traits::{bool#8}]
+ Source: 'src/traits.rs', lines 174:0-174:29 -/
def traits.WithConstTyBool32Inst : WithConstTy Bool 32#usize := {
LEN1 := bool_len1_c
LEN2 := with_const_ty_len2_c
@@ -232,153 +275,183 @@ def traits.WithConstTyBool32Inst : WithConstTy Bool 32#usize := {
f := Bool.f
}
-/- [traits::use_with_const_ty1]: forward function -/
+/- [traits::use_with_const_ty1]: forward function
+ Source: 'src/traits.rs', lines 183:0-183:75 -/
def use_with_const_ty1
(H : Type) (LEN : Usize) (inst : WithConstTy H LEN) : Result Usize :=
let i := inst.LEN1
Result.ret i
-/- [traits::use_with_const_ty2]: forward function -/
+/- [traits::use_with_const_ty2]: forward function
+ Source: 'src/traits.rs', lines 187:0-187:73 -/
def use_with_const_ty2
(H : Type) (LEN : Usize) (inst : WithConstTy H LEN) (w : inst.W) :
Result Unit
:=
Result.ret ()
-/- [traits::use_with_const_ty3]: forward function -/
+/- [traits::use_with_const_ty3]: forward function
+ Source: 'src/traits.rs', lines 189:0-189:80 -/
def use_with_const_ty3
(H : Type) (LEN : Usize) (inst : WithConstTy H LEN) (x : inst.W) :
Result U64
:=
inst.W_clause_0.to_u64 x
-/- [traits::test_where1]: forward function -/
+/- [traits::test_where1]: forward function
+ Source: 'src/traits.rs', lines 193:0-193:40 -/
def test_where1 (T : Type) (_x : T) : Result Unit :=
Result.ret ()
-/- [traits::test_where2]: forward function -/
+/- [traits::test_where2]: forward function
+ Source: 'src/traits.rs', lines 194:0-194:57 -/
def test_where2
(T : Type) (inst : WithConstTy T 32#usize) (_x : U32) : Result Unit :=
Result.ret ()
-/- [alloc::string::String] -/
+/- [alloc::string::String]
+ Source: '/rustc/d59363ad0b6391b7fc5bbb02c9ccf9300eef3753/library/alloc/src/string.rs', lines 365:0-365:17 -/
axiom alloc.string.String : Type
-/- Trait declaration: [traits::ParentTrait0] -/
+/- Trait declaration: [traits::ParentTrait0]
+ Source: 'src/traits.rs', lines 200:0-200:22 -/
structure ParentTrait0 (Self : Type) where
W : Type
get_name : Self → Result alloc.string.String
get_w : Self → Result W
-/- Trait declaration: [traits::ParentTrait1] -/
+/- Trait declaration: [traits::ParentTrait1]
+ Source: 'src/traits.rs', lines 205:0-205:22 -/
structure ParentTrait1 (Self : Type) where
-/- Trait declaration: [traits::ChildTrait] -/
+/- Trait declaration: [traits::ChildTrait]
+ Source: 'src/traits.rs', lines 206:0-206:49 -/
structure ChildTrait (Self : Type) where
parent_clause_0 : ParentTrait0 Self
parent_clause_1 : ParentTrait1 Self
-/- [traits::test_child_trait1]: forward function -/
+/- [traits::test_child_trait1]: forward function
+ Source: 'src/traits.rs', lines 209:0-209:56 -/
def test_child_trait1
(T : Type) (inst : ChildTrait T) (x : T) : Result alloc.string.String :=
inst.parent_clause_0.get_name x
-/- [traits::test_child_trait2]: forward function -/
+/- [traits::test_child_trait2]: forward function
+ Source: 'src/traits.rs', lines 213:0-213:54 -/
def test_child_trait2
(T : Type) (inst : ChildTrait T) (x : T) : Result inst.parent_clause_0.W :=
inst.parent_clause_0.get_w x
-/- [traits::order1]: forward function -/
+/- [traits::order1]: forward function
+ Source: 'src/traits.rs', lines 219:0-219:59 -/
def order1
(T U : Type) (inst : ParentTrait0 T) (inst0 : ParentTrait0 U) :
Result Unit
:=
Result.ret ()
-/- Trait declaration: [traits::ChildTrait1] -/
+/- Trait declaration: [traits::ChildTrait1]
+ Source: 'src/traits.rs', lines 222:0-222:35 -/
structure ChildTrait1 (Self : Type) where
parent_clause_0 : ParentTrait1 Self
-/- Trait implementation: [traits::{usize#9}] -/
+/- Trait implementation: [traits::{usize#9}]
+ Source: 'src/traits.rs', lines 224:0-224:27 -/
def traits.ParentTrait1UsizeInst : ParentTrait1 Usize := {
}
-/- Trait implementation: [traits::{usize#10}] -/
+/- Trait implementation: [traits::{usize#10}]
+ Source: 'src/traits.rs', lines 225:0-225:26 -/
def traits.ChildTrait1UsizeInst : ChildTrait1 Usize := {
parent_clause_0 := traits.ParentTrait1UsizeInst
}
-/- Trait declaration: [traits::Iterator] -/
+/- Trait declaration: [traits::Iterator]
+ Source: 'src/traits.rs', lines 229:0-229:18 -/
structure Iterator (Self : Type) where
Item : Type
-/- Trait declaration: [traits::IntoIterator] -/
+/- Trait declaration: [traits::IntoIterator]
+ Source: 'src/traits.rs', lines 233:0-233:22 -/
structure IntoIterator (Self : Type) where
Item : Type
IntoIter : Type
IntoIter_clause_0 : Iterator IntoIter
into_iter : Self → Result IntoIter
-/- Trait declaration: [traits::FromResidual] -/
+/- Trait declaration: [traits::FromResidual]
+ Source: 'src/traits.rs', lines 250:0-250:21 -/
structure FromResidual (Self T : Type) where
-/- Trait declaration: [traits::Try] -/
+/- Trait declaration: [traits::Try]
+ Source: 'src/traits.rs', lines 246:0-246:48 -/
structure Try (Self : Type) where
Residual : Type
parent_clause_0 : FromResidual Self Residual
-/- Trait declaration: [traits::WithTarget] -/
+/- Trait declaration: [traits::WithTarget]
+ Source: 'src/traits.rs', lines 252:0-252:20 -/
structure WithTarget (Self : Type) where
Target : Type
-/- Trait declaration: [traits::ParentTrait2] -/
+/- Trait declaration: [traits::ParentTrait2]
+ Source: 'src/traits.rs', lines 256:0-256:22 -/
structure ParentTrait2 (Self : Type) where
U : Type
U_clause_0 : WithTarget U
-/- Trait declaration: [traits::ChildTrait2] -/
+/- Trait declaration: [traits::ChildTrait2]
+ Source: 'src/traits.rs', lines 260:0-260:35 -/
structure ChildTrait2 (Self : Type) where
parent_clause_0 : ParentTrait2 Self
convert : parent_clause_0.U → Result parent_clause_0.U_clause_0.Target
-/- Trait implementation: [traits::{u32#11}] -/
+/- Trait implementation: [traits::{u32#11}]
+ Source: 'src/traits.rs', lines 264:0-264:23 -/
def traits.WithTargetU32Inst : WithTarget U32 := {
Target := U32
}
-/- Trait implementation: [traits::{u32#12}] -/
+/- Trait implementation: [traits::{u32#12}]
+ Source: 'src/traits.rs', lines 268:0-268:25 -/
def traits.ParentTrait2U32Inst : ParentTrait2 U32 := {
U := U32
U_clause_0 := traits.WithTargetU32Inst
}
-/- [traits::{u32#13}::convert]: forward function -/
+/- [traits::{u32#13}::convert]: forward function
+ Source: 'src/traits.rs', lines 273:4-273:29 -/
def U32.convert (x : U32) : Result U32 :=
Result.ret x
-/- Trait implementation: [traits::{u32#13}] -/
+/- Trait implementation: [traits::{u32#13}]
+ Source: 'src/traits.rs', lines 272:0-272:24 -/
def traits.ChildTrait2U32Inst : ChildTrait2 U32 := {
parent_clause_0 := traits.ParentTrait2U32Inst
convert := U32.convert
}
-/- Trait declaration: [traits::CFnOnce] -/
+/- Trait declaration: [traits::CFnOnce]
+ Source: 'src/traits.rs', lines 286:0-286:23 -/
structure CFnOnce (Self Args : Type) where
Output : Type
call_once : Self → Args → Result Output
-/- Trait declaration: [traits::CFnMut] -/
+/- Trait declaration: [traits::CFnMut]
+ Source: 'src/traits.rs', lines 292:0-292:37 -/
structure CFnMut (Self Args : Type) where
parent_clause_0 : CFnOnce Self Args
call_mut : Self → Args → Result parent_clause_0.Output
call_mut_back : Self → Args → parent_clause_0.Output → Result Self
-/- Trait declaration: [traits::CFn] -/
+/- Trait declaration: [traits::CFn]
+ Source: 'src/traits.rs', lines 296:0-296:33 -/
structure CFn (Self Args : Type) where
parent_clause_0 : CFnMut Self Args
call_mut : Self → Args → Result parent_clause_0.parent_clause_0.Output
-/- [traits::incr_u32]: forward function -/
+/- [traits::incr_u32]: forward function
+ Source: 'src/traits.rs', lines 300:0-300:30 -/
def incr_u32 (x : U32) : Result U32 :=
x + 1#u32