File tree Expand file tree Collapse file tree 1 file changed +34
-0
lines changed
Expand file tree Collapse file tree 1 file changed +34
-0
lines changed Original file line number Diff line number Diff line change 1+ example (n : Nat)
2+ (f : Nat → Rat → Rat)
3+ (x : Rat)
4+ (H : ∀ (x : Rat), 0 ≤ x →
5+ (4 < x → f n x < 2 * x) ∧ (x = 4 → f n x = 2 * x) ∧ (x < 4 → 2 * x < f n x)) :
6+ x ∈ [4 ] ↔ f n x = 2 * x := by
7+ fail_if_success grind
8+ sorry
9+
10+ example (n : Nat)
11+ (f : Nat → Rat → Rat)
12+ (x : Rat)
13+ (_ : x ≥ 0 )
14+ (H : ∀ (x : Rat), 0 ≤ x →
15+ (4 < x → f n x < 2 * x) ∧ (x = 4 → f n x = 2 * x) ∧ (x < 4 → 2 * x < f n x)) :
16+ x ∈ [4 ] ↔ f n x = 2 * x := by
17+ grind
18+
19+ example (n : Nat)
20+ (f : Nat → Rat → Rat)
21+ (x : Rat)
22+ (_ : x ≥ 0 )
23+ (H : ∀ (x : Rat), 0 ≤ x →
24+ (4 < x → f n x < 2 * x) ∧ (x = 4 → f n x = 2 * x) ∧ (x < 4 → 2 * x < f n x)) :
25+ f n x = 2 * x → x ∈ [4 ] := by
26+ grind
27+
28+ example (n : Nat)
29+ (f : Nat → Rat → Rat)
30+ (x : Rat)
31+ (H : ∀ (x : Rat), 0 ≤ x →
32+ (4 < x → f n x < 2 * x) ∧ (x = 4 → f n x = 2 * x) ∧ (x < 4 → 2 * x < f n x)) :
33+ x ∈ [4 ] → f n x = 2 * x := by
34+ grind
You can’t perform that action at this time.
0 commit comments