File tree Expand file tree Collapse file tree 1 file changed +15
-0
lines changed Expand file tree Collapse file tree 1 file changed +15
-0
lines changed Original file line number Diff line number Diff line change @@ -70,6 +70,21 @@ testIndep 6 50 by
70
70
trivial
71
71
-/
72
72
73
+ /--
74
+ #### Independent rules.
75
+
76
+ This test compares the efficiency of the procedures on independent rules
77
+ and hypotheses.
78
+
79
+ Consider a set of propositions `P := {Pᵢⱼ | 1 ≤ i ≤ nRs and 1 ≤ j ≤ nPs}` and
80
+ `Q := {Qᵢ | 1 ≤ i ≤ nRs}`.
81
+ We run the procedures we with the `nRs` following rules `rᵢ : Pᵢ₁ → ... → Pᵢₙₚₛ → Qᵢ`
82
+ and a context containing precisely `P`.
83
+
84
+ - `nPs` : Number of premises in the rules.
85
+ - `nRs` : Number of unique rules; they are independent but have the same number
86
+ of premises.
87
+ -/
73
88
def runTestIndep (nPs : Nat) (nRs : Nat) : CommandElabM Nanos := do
74
89
let mut nPs := Syntax.mkNatLit nPs
75
90
let mut nRs := Syntax.mkNatLit nRs
You can’t perform that action at this time.
0 commit comments