diff -r 50d3059de9c6 -r 6e2479089226 ProgTutorial/Base.thy --- a/ProgTutorial/Base.thy Tue May 14 13:39:31 2019 +0200 +++ b/ProgTutorial/Base.thy Tue May 14 16:59:53 2019 +0200 @@ -3,17 +3,12 @@ "~~/src/HOL/Library/LaTeXsugar" begin -ML \@{assert} true\ -ML \@{print} (2 + 3 +4)\ - +print_ML_antiquotations -print_ML_antiquotations -text \ -Can we put an ML-val into the text? +text \Hallo ML Antiquotation: +@{ML \2 + 3\} +\ -@{ML [display] \2 + 3\} - -\ notation (latex output) Cons ("_ # _" [66,65] 65) @@ -30,17 +25,16 @@ HOLogic.mk_Trueprop (HOLogic.mk_imp (lhs n n, rhs n))*} ML_file "output_tutorial.ML" -text \ -Can we put an ML-val into the text? - -@{ML [gray] \2 + 3\} -\ - ML_file "antiquote_setup.ML" (*setup {* OutputTutorial.setup *}*) (* Seems to be standard now, we don't need this anymoe *) setup {* AntiquoteSetup.setup *} +print_ML_antiquotations + +text \Hallo ML Antiquotation: +@{ML \2 + 3\ } +\ end \ No newline at end of file