doc-src/IsarImplementation/Thy/Base.thy
author wenzelm
Thu, 21 Oct 2010 20:00:46 +0100
changeset 39876 1ff9bce085bd
parent 39866 5ec01d5acd0c
child 40110 93e7935d4cb5
permissions -rw-r--r--
preliminary material on "Concrete syntax and type-checking";

theory Base
imports Main
uses "../../antiquote_setup.ML"
begin

(* FIXME move to src/Pure/ML/ml_antiquote.ML *)
ML {*
  ML_Antiquote.inline "assert"
    (Scan.succeed "(fn b => if b then () else raise General.Fail \"Assertion failed\")")
*}

end