author | Norbert Schirmer <norbert.schirmer@web.de> |
Wed, 22 May 2019 13:24:30 +0200 | |
changeset 575 | c3dbc04471a9 |
parent 573 | 321e220a6baa |
permissions | -rw-r--r-- |
23 | 1 |
theory Base |
459 | 2 |
imports Main |
3 |
"~~/src/HOL/Library/LaTeXsugar" |
|
23 | 4 |
begin |
5 |
||
573
321e220a6baa
accomodate to upcoming Isabelle 2019
Norbert Schirmer <norbert.schirmer@web.de>
parents:
572
diff
changeset
|
6 |
|
394 | 7 |
notation (latex output) |
8 |
Cons ("_ # _" [66,65] 65) |
|
9 |
||
565
cecd7a941885
isabelle update_cartouches -t
Norbert Schirmer <norbert.schirmer@web.de>
parents:
564
diff
changeset
|
10 |
ML %linenosgrayML\<open>fun P n = @{term "P::nat \<Rightarrow> bool"} $ (HOLogic.mk_number @{typ "nat"} n) |
396 | 11 |
|
12 |
fun rhs 1 = P 1 |
|
13 |
| rhs n = HOLogic.mk_conj (P n, rhs (n - 1)) |
|
14 |
||
15 |
fun lhs 1 n = HOLogic.mk_imp (HOLogic.mk_eq (P 1, P n), rhs n) |
|
16 |
| lhs m n = HOLogic.mk_conj (HOLogic.mk_imp |
|
17 |
(HOLogic.mk_eq (P (m - 1), P m), rhs n), lhs (m - 1) n) |
|
18 |
||
19 |
fun de_bruijn n = |
|
565
cecd7a941885
isabelle update_cartouches -t
Norbert Schirmer <norbert.schirmer@web.de>
parents:
564
diff
changeset
|
20 |
HOLogic.mk_Trueprop (HOLogic.mk_imp (lhs n n, rhs n))\<close> |
346
0fea8b7a14a1
tuned the ML-output mechanism; tuned slightly the text
Christian Urban <urbanc@in.tum.de>
parents:
328
diff
changeset
|
21 |
|
538
e9fd5eff62c1
removed "use" for "ML_file"
Christian Urban <urbanc@in.tum.de>
parents:
535
diff
changeset
|
22 |
ML_file "output_tutorial.ML" |
e9fd5eff62c1
removed "use" for "ML_file"
Christian Urban <urbanc@in.tum.de>
parents:
535
diff
changeset
|
23 |
ML_file "antiquote_setup.ML" |
346
0fea8b7a14a1
tuned the ML-output mechanism; tuned slightly the text
Christian Urban <urbanc@in.tum.de>
parents:
328
diff
changeset
|
24 |
|
565
cecd7a941885
isabelle update_cartouches -t
Norbert Schirmer <norbert.schirmer@web.de>
parents:
564
diff
changeset
|
25 |
setup \<open>AntiquoteSetup.setup\<close> |
346
0fea8b7a14a1
tuned the ML-output mechanism; tuned slightly the text
Christian Urban <urbanc@in.tum.de>
parents:
328
diff
changeset
|
26 |
|
239
b63c72776f03
replaced "warning" with "writeln"
Christian Urban <urbanc@in.tum.de>
parents:
224
diff
changeset
|
27 |
end |